src/HOL/W0/Maybe.ML
changeset 4831 dae4d63a1318
parent 4089 96fba19bcbe2
child 5069 3ea049f7979d
--- a/src/HOL/W0/Maybe.ML	Mon Apr 27 16:45:11 1998 +0200
+++ b/src/HOL/W0/Maybe.ML	Mon Apr 27 16:45:27 1998 +0200
@@ -16,17 +16,17 @@
 
 Addsimps [bind_Ok,bind_Fail];
 
-(* expansion of bind *)
+(* case splitting of bind *)
 goal thy
   "P(res bind f) = ((res = Fail --> P Fail) & (!s. res = Ok s --> P(f s)))";
-by (maybe.induct_tac "res" 1);
+by (induct_tac "res" 1);
 by (fast_tac (HOL_cs addss simpset()) 1);
 by (Asm_simp_tac 1);
-qed "expand_bind";
+qed "split_bind";
 
 goal Maybe.thy
   "((m bind f) = Fail) = ((m=Fail) | (? p. m = Ok p & f p = Fail))";
-by (simp_tac (simpset() addsplits [expand_bind]) 1);
+by (simp_tac (simpset() addsplits [split_bind]) 1);
 qed "bind_eq_Fail";
 
 Addsimps [bind_eq_Fail];