diff -r 56057198e4f5 -r 70c10dc41606 thys3/FBound.thy --- a/thys3/FBound.thy Fri May 26 08:09:30 2023 +0100 +++ b/thys3/FBound.thy Fri May 26 08:10:17 2023 +0100 @@ -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)"