test/Tools/isac/Test_Theory.thy
author wneuper <Walther.Neuper@jku.at>
Wed, 27 Sep 2023 12:17:44 +0200
changeset 60755 b817019bfda7
parent 60753 30eb1f314f5c
child 60760 3b173806efe2
permissions -rw-r--r--
prepare 9: I_Model.complete* all replaced by I_Model.s_make_complete
wneuper@59119
     1
(* use this theory for tests before Build_Isac.thy has succeeded *)
Walther@60576
     2
theory Test_Theory imports "$ISABELLE_ISAC/Build_Isac"
Walther@60736
     3
  "$ISABELLE_ISAC_TEST/Tools/isac/Specify/refine"        (* setup for refine.sml   *)
neuper@52102
     4
begin                                                                            
wenzelm@60192
     5
ML_file "$ISABELLE_ISAC/BaseDefinitions/libraryC.sml"
neuper@52102
     6
wneuper@59472
     7
section \<open>code for copy & paste ===============================================================\<close>
Walther@60737
     8
text \<open>
Walther@60737
     9
  declare [[show_types]] 
Walther@60737
    10
  declare [[show_sorts]]
Walther@60737
    11
  find_theorems "?a <= ?a"
Walther@60737
    12
  
Walther@60737
    13
  print_theorems
Walther@60737
    14
  print_facts
Walther@60737
    15
  print_statement ""
Walther@60737
    16
  print_theory
Walther@60737
    17
  ML_command \<open>Pretty.writeln prt\<close>
Walther@60737
    18
  declare [[ML_print_depth = 999]]
Walther@60737
    19
  declare [[ML_exception_trace]]
Walther@60737
    20
\<close>
Walther@60751
    21
(** )
Walther@60751
    22
  (@{print} {a = "dict_cond_ord ([], [])"}; EQUAL)
Walther@60751
    23
( **)
wneuper@59472
    24
ML \<open>
Walther@60710
    25
\<close> ML \<open>
walther@59686
    26
"~~~~~ fun xxx , args:"; val () = ();
walther@59686
    27
"~~~~~ and xxx , args:"; val () = ();
Walther@60576
    28
"~~~~~ from fun xxx \<longrightarrow>fun yyy \<longrightarrow>fun zzz , return:"; val () = ();
Walther@60576
    29
"~~~~~ continue fun xxx"; val () = ();
Walther@60729
    30
(*if*) (*then*); (*else*); (*andalso*)  (*case*) (*of*);  (*return value*); (*in*) (*end*);
walther@59686
    31
"xx"
Walther@60629
    32
^ "xxx"   (*+*) (*+++*) (*keep for continuing YYYYY*) (*isa*) (*isa2*) (**)
Walther@60729
    33
\<close> ML \<open> (*//----------- build fun XXXXX -----------------------------------------------------\\*)
Walther@60729
    34
(*//------------------ build fun XXXXX -----------------------------------------------------\\*)
Walther@60729
    35
(*\\------------------ build fun XXXXX -----------------------------------------------------//*)
Walther@60729
    36
\<close> ML \<open> (*\\----------- build fun XXXXX -----------------------------------------------------//*)
Walther@60737
    37
Walther@60751
    38
\<close> ML \<open> (*//----------- setup test data for XXXXX -------------------------------------------\\*)
Walther@60751
    39
(*//------------------ setup test data for XXXXX -------------------------------------------\\*)
Walther@60751
    40
(*\\------------------ setup test data for XXXXX -------------------------------------------//*)
Walther@60751
    41
\<close> ML \<open> (*\\----------- setup test data for XXXXX -------------------------------------------//*)
Walther@60751
    42
Walther@60682
    43
val return_XXXXX = "XXXXX"
Walther@60576
    44
\<close> ML \<open> (*//----------- step into XXXXX -----------------------------------------------------\\*)
Walther@60576
    45
(*//------------------ step into XXXXX -----------------------------------------------------\\*)
Walther@60715
    46
\<close> ML \<open> (*||----------- contine XXXXX ---------------------------------------------------------*)
Walther@60715
    47
(*||------------------ contine XXXXX ---------------------------------------------------------*)
Walther@60576
    48
(*\\------------------ step into XXXXX -----------------------------------------------------//*)
Walther@60576
    49
\<close> ML \<open> (*\\----------- step into XXXXX -----------------------------------------------------//*)
Walther@60710
    50
val "XXXXX" = return_XXXXX;
Walther@60576
    51
Walther@60576
    52
(* final test ... ----------------------------------------------------------------------------*)
Walther@60576
    53
Walther@60576
    54
\<close> ML \<open> (*//----------- inserted hidden code ------------------------------------------------\\*)
Walther@60576
    55
(*//------------------ inserted hidden code ------------------------------------------------\\*)
Walther@60576
    56
(*\\------------------ inserted hidden code ------------------------------------------------//*)
Walther@60576
    57
\<close> ML \<open> (*\\----------- inserted hidden code ------------------------------------------------//*)
Walther@60576
    58
walther@59723
    59
\<close> ML \<open>
wneuper@59472
    60
\<close>
neuper@52102
    61
Walther@60658
    62
section \<open>===================================================================================\<close>
Walther@60725
    63
section \<open>=====  ============================================================================\<close>
wneuper@59472
    64
ML \<open>
wneuper@59472
    65
\<close> ML \<open>
Walther@60733
    66
Walther@60733
    67
\<close> ML \<open>
Walther@60733
    68
\<close>
Walther@60733
    69
Walther@60733
    70
section \<open>===================================================================================\<close>
Walther@60755
    71
section \<open>=====  ============================================================================\<close>
Walther@60733
    72
ML \<open>
Walther@60736
    73
\<close> ML \<open>
Walther@60752
    74
Walther@60752
    75
\<close> ML \<open>
Walther@60752
    76
\<close>
Walther@60752
    77
Walther@60752
    78
section \<open>===================================================================================\<close>
Walther@60736
    79
section \<open>=====   ===========================================================================\<close>
Walther@60736
    80
ML \<open>
Walther@60715
    81
\<close> ML \<open>
Walther@60715
    82
Walther@60723
    83
\<close> ML \<open>
Walther@60736
    84
\<close>
Walther@60736
    85
neuper@52102
    86
end