We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent f87573d commit f6a7e00Copy full SHA for f6a7e00
src/coalgebras/itreeTauScript.sml
@@ -1166,11 +1166,11 @@ QED
1166
(* coinduction upto stripping finite taus, useful for iter and friends *)
1167
Inductive after_taus:
1168
[~rel:]
1169
- (R x y ==> after_taus R x y) /\
+ (R x y ==> after_taus R x y)
1170
[~tauL:]
1171
- (after_taus R x y ==> after_taus R (Tau x) y) /\
+ (after_taus R x y ==> after_taus R (Tau x) y)
1172
[~tauR:]
1173
- (after_taus R x y ==> after_taus R x (Tau y)) /\
+ (after_taus R x y ==> after_taus R x (Tau y))
1174
[~vis:]
1175
((!r. after_taus R (k r) (k' r)) ==> after_taus R (Vis e k) (Vis e k'))
1176
End
0 commit comments