| author | blanchet | 
| Thu, 05 May 2011 12:40:48 +0200 | |
| changeset 42699 | d4f5fec71ded | 
| parent 41959 | b460124855b8 | 
| permissions | -rw-r--r-- | 
| 41959 | 1 | (* Title: HOL/Matrix/Compute_Oracle/Compute_Oracle.thy | 
| 23173 
51179ca0c429
proper theory setup for compute oracle (based on CPure);
 wenzelm parents: diff
changeset | 2 | Author: Steven Obua, TU Munich | 
| 
51179ca0c429
proper theory setup for compute oracle (based on CPure);
 wenzelm parents: diff
changeset | 3 | |
| 
51179ca0c429
proper theory setup for compute oracle (based on CPure);
 wenzelm parents: diff
changeset | 4 | Steven Obua's evaluator. | 
| 
51179ca0c429
proper theory setup for compute oracle (based on CPure);
 wenzelm parents: diff
changeset | 5 | *) | 
| 
51179ca0c429
proper theory setup for compute oracle (based on CPure);
 wenzelm parents: diff
changeset | 6 | |
| 37869 | 7 | theory Compute_Oracle imports HOL | 
| 25217 | 8 | uses "am.ML" "am_compiler.ML" "am_interpreter.ML" "am_ghc.ML" "am_sml.ML" "report.ML" "compute.ML" "linker.ML" | 
| 23173 
51179ca0c429
proper theory setup for compute oracle (based on CPure);
 wenzelm parents: diff
changeset | 9 | begin | 
| 
51179ca0c429
proper theory setup for compute oracle (based on CPure);
 wenzelm parents: diff
changeset | 10 | |
| 23663 | 11 | end |