diff -r cf7a5c863831 -r 6c13f76c070b thys3/FBound.thy --- a/thys3/FBound.thy Wed Feb 15 11:52:22 2023 +0000 +++ b/thys3/FBound.thy Thu Feb 16 23:23:22 2023 +0000 @@ -18,6 +18,7 @@ | "rerase (AALTs bs rs) = RALTS (map rerase rs)" | "rerase (ASEQ _ r1 r2) = RSEQ (rerase r1) (rerase r2)" | "rerase (ASTAR _ r) = RSTAR (rerase r)" +| "rerase (ANTIMES _ r n) = RNTIMES (rerase r) n" lemma eq1_rerase: shows "x ~1 y \ (rerase x) = (rerase y)"