| author | paulson | 
| Mon, 24 May 1999 15:53:28 +0200 | |
| changeset 6715 | 89891b0b596f | 
| parent 6466 | 2eba94dc5951 | 
| child 7295 | fe09a0c5cebe | 
| permissions | -rw-r--r-- | 
(* Title: HOL/Modelcheck/MuckeExample2.ML ID: $Id$ Author: Olaf Mueller, Jan Philipps, Robert Sandner Copyright 1997 TU Muenchen *) (* prints the mucke output on the screen *) (* trace_mc := true; *) val Reach_rws = [Init_def,R_def,Reach_def,Reach2_def]; (* goal thy "Reach2 True"; by (simp_tac (Mucke_ss addsimps Reach_rws) 1); by (mc_mucke_tac thy [] 1); qed "Reach_thm"; (* Alternative: *) goal thy "Reach2 True"; by (mc_mucke_tac thy Reach_rws 1); qed "Reach_thm"; *)